# HG changeset patch # User Cezary Kaliszyk # Date 1264677889 -3600 # Node ID 9d35c6145dd208f9123609209a477b6762fabaec # Parent a88e16b69d0f891143f32579e7b0581aa30f45c2 Renamed Bexeq to Bex1_rel diff -r a88e16b69d0f -r 9d35c6145dd2 Attic/Unused.thy --- a/Attic/Unused.thy Thu Jan 28 10:52:10 2010 +0100 +++ b/Attic/Unused.thy Thu Jan 28 12:24:49 2010 +0100 @@ -6,9 +6,9 @@ by(auto simp add: QUOT_TRUE_def) syntax - "Bexeq" :: "id \ ('a \ 'a \ bool) \ ('a \ bool) \ bool" ("(3\!!_\_./ _)" [0, 0, 10] 10) + "Bex1_rel" :: "id \ ('a \ 'a \ bool) \ ('a \ bool) \ bool" ("(3\!!_\_./ _)" [0, 0, 10] 10) translations - "\!!x\A. P" == "Bexeq A (%x. P)" + "\!!x\A. P" == "Bex1_rel A (%x. P)" (* Atomize infrastructure *) diff -r a88e16b69d0f -r 9d35c6145dd2 Quot/Examples/SigmaEx.thy --- a/Quot/Examples/SigmaEx.thy Thu Jan 28 10:52:10 2010 +0100 +++ b/Quot/Examples/SigmaEx.thy Thu Jan 28 12:24:49 2010 +0100 @@ -128,8 +128,8 @@ sorry -lemma bex1_bex1reg: "(\!x\Respects R. P x) \ (Bexeq R (\x. P x))" -apply (simp add: Bex1_def Ex1_def Bexeq_def in_respects) +lemma bex1_bex1reg: "(\!x\Respects R. P x) \ (Bex1_rel R (\x. P x))" +apply (simp add: Bex1_def Ex1_def Bex1_rel_def in_respects) apply clarify apply auto apply (rule bexI) @@ -207,10 +207,10 @@ \ fpar\Respects (op = ===> op = ===> alpha_method ===> op =). \ fsgm\Respects (op = ===> (op = ===> alpha_obj) ===> op =). - Bexeq (alpha_obj ===> op =) (\hom_o\robj \ 'a . - Bexeq (list_rel (prod_rel (op =) alpha_method) ===> op =) (\hom_d\(char list \ rmethod) list \ 'b. - Bexeq ((prod_rel (op =) alpha_method) ===> op =) (\hom_e\char list \ rmethod \ 'c. - Bexeq (alpha_method ===> op =) (\hom_m\rmethod \ 'd. + Bex1_rel (alpha_obj ===> op =) (\hom_o\robj \ 'a . + Bex1_rel (list_rel (prod_rel (op =) alpha_method) ===> op =) (\hom_d\(char list \ rmethod) list \ 'b. + Bex1_rel ((prod_rel (op =) alpha_method) ===> op =) (\hom_e\char list \ rmethod \ 'c. + Bex1_rel (alpha_method ===> op =) (\hom_m\rmethod \ 'd. ( (\x. hom_o (rVar x) = fvar x) \ (\d. hom_o (rObj d) = fobj (hom_d d) d) \ diff -r a88e16b69d0f -r 9d35c6145dd2 Quot/QuotBase.thy --- a/Quot/QuotBase.thy Thu Jan 28 10:52:10 2010 +0100 +++ b/Quot/QuotBase.thy Thu Jan 28 12:24:49 2010 +0100 @@ -451,19 +451,19 @@ using a unfolding Quotient_def Bex_def in_respects fun_map_def id_apply by metis -section {* Bexeq quantifier *} +section {* Bex1_rel quantifier *} definition - Bexeq :: "('a \ 'a \ bool) \ ('a \ bool) \ bool" + Bex1_rel :: "('a \ 'a \ bool) \ ('a \ bool) \ bool" where - "Bexeq R P \ (\x \ Respects R. P x) \ (\x \ Respects R. \y \ Respects R. ((P x \ P y) \ (R x y)))" + "Bex1_rel R P \ (\x \ Respects R. P x) \ (\x \ Respects R. \y \ Respects R. ((P x \ P y) \ (R x y)))" (* TODO/FIXME: simplify the repetitions in this proof *) lemma bexeq_rsp: assumes a: "Quotient R absf repf" - shows "((R ===> op =) ===> op =) (Bexeq R) (Bexeq R)" + shows "((R ===> op =) ===> op =) (Bex1_rel R) (Bex1_rel R)" apply simp -unfolding Bexeq_def +unfolding Bex1_rel_def apply rule apply rule apply rule @@ -500,9 +500,9 @@ lemma ex1_prs: assumes a: "Quotient R absf repf" - shows "((absf ---> id) ---> id) (Bexeq R) f = Ex1 f" + shows "((absf ---> id) ---> id) (Bex1_rel R) f = Ex1 f" apply simp -apply (subst Bexeq_def) +apply (subst Bex1_rel_def) apply (subst Bex_def) apply (subst Ex1_def) apply simp @@ -535,8 +535,8 @@ apply metis done -lemma bex1_bexeq_reg: "(\!x\Respects R. P x) \ (Bexeq R (\x. P x))" - apply (simp add: Bex1_def Ex1_def Bexeq_def in_respects) +lemma bex1_bexeq_reg: "(\!x\Respects R. P x) \ (Bex1_rel R (\x. P x))" + apply (simp add: Bex1_def Ex1_def Bex1_rel_def in_respects) apply clarify apply auto apply (rule bexI) diff -r a88e16b69d0f -r 9d35c6145dd2 Quot/quotient_tacs.ML --- a/Quot/quotient_tacs.ML Thu Jan 28 10:52:10 2010 +0100 +++ b/Quot/quotient_tacs.ML Thu Jan 28 12:24:49 2010 +0100 @@ -366,7 +366,7 @@ => rtac @{thm fun_rel_id} THEN' quot_true_tac ctxt unlam | (Const (@{const_name fun_rel}, _) $ _ $ _) $ - (Const(@{const_name Bexeq},_) $ _) $ (Const(@{const_name Bexeq},_) $ _) + (Const(@{const_name Bex1_rel},_) $ _) $ (Const(@{const_name Bex1_rel},_) $ _) => rtac @{thm bexeq_rsp} THEN' quotient_tac ctxt | (_ $