Skip to content
Snippets Groups Projects
Commit 9af65178 authored by Robbert Krebbers's avatar Robbert Krebbers
Browse files

Make Program obligations Transparent by default.

This may save the need to seal off some stuff.
parent 8759beb5
No related branches found
No related tags found
No related merge requests found
...@@ -148,8 +148,8 @@ Arguments agreeC : clear implicits. ...@@ -148,8 +148,8 @@ Arguments agreeC : clear implicits.
Arguments agreeR : clear implicits. Arguments agreeR : clear implicits.
Program Definition agree_map {A B} (f : A B) (x : agree A) : agree B := Program Definition agree_map {A B} (f : A B) (x : agree A) : agree B :=
{| agree_car n := f (x n); agree_is_valid := agree_is_valid x |}. {| agree_car n := f (x n); agree_is_valid := agree_is_valid x;
Solve Obligations with auto using agree_valid_S. agree_valid_S := agree_valid_S _ x |}.
Lemma agree_map_id {A} (x : agree A) : agree_map id x = x. Lemma agree_map_id {A} (x : agree A) : agree_map id x = x.
Proof. by destruct x. Qed. Proof. by destruct x. Qed.
Lemma agree_map_compose {A B C} (f : A B) (g : B C) (x : agree A) : Lemma agree_map_compose {A B C} (f : A B) (g : B C) (x : agree A) :
......
...@@ -7,6 +7,7 @@ structures. *) ...@@ -7,6 +7,7 @@ structures. *)
Global Generalizable All Variables. Global Generalizable All Variables.
Global Set Automatic Coercions Import. Global Set Automatic Coercions Import.
Global Set Asymmetric Patterns. Global Set Asymmetric Patterns.
Global Unset Transparent Obligations.
From Coq Require Export Morphisms RelationClasses List Bool Utf8 Program Setoid. From Coq Require Export Morphisms RelationClasses List Bool Utf8 Program Setoid.
Obligation Tactic := idtac. Obligation Tactic := idtac.
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment