Normalise equation only for morphism, not thm stored in theory.
authorballarin
Sun, 29 Mar 2009 17:22:17 +0200
changeset 30781 7fb900cad123
parent 30780 c3f1e8a9e0b5
child 30782 38e477e8524f
Normalise equation only for morphism, not thm stored in theory.
src/Pure/Isar/expression.ML
--- a/src/Pure/Isar/expression.ML	Sat Mar 28 22:14:21 2009 +0100
+++ b/src/Pure/Isar/expression.ML	Sun Mar 29 17:22:17 2009 +0200
@@ -833,10 +833,10 @@
                Locale.activate_global_facts (name, morph $> export)) regs
       | store_eqns_activate regs eqs thy =
           let
-            val eqs' = eqs |> map (Morphism.thm (export' $> export) #>
-              LocalDefs.meta_rewrite_rule (ProofContext.init thy) #>
+            val eqs' = eqs |> map (Morphism.thm (export' $> export));
+            val morph_eqs = eqs' |> map (LocalDefs.meta_rewrite_rule (ProofContext.init thy) #>
               Drule.abs_def);
-            val eq_morph = Element.eq_morphism thy eqs';
+            val eq_morph = Element.eq_morphism thy morph_eqs;
             val eq_attns' = map ((apsnd o map) (Attrib.attribute_i thy)) eq_attns;
           in
             thy