src/ZF/Datatype_ZF.thy
changeset 51930 52fd62618631
parent 51717 9e7d1c139569
child 54388 8b165615ffe3
--- a/src/ZF/Datatype_ZF.thy	Sat May 11 16:13:08 2013 +0200
+++ b/src/ZF/Datatype_ZF.thy	Sat May 11 16:57:18 2013 +0200
@@ -81,9 +81,9 @@
        val lname = #1 (dest_Const lhead) handle TERM _ => raise Match;
        val rname = #1 (dest_Const rhead) handle TERM _ => raise Match;
        val lcon_info = the (Symtab.lookup (ConstructorsData.get thy) lname)
-         handle Option => raise Match;
+         handle Option.Option => raise Match;
        val rcon_info = the (Symtab.lookup (ConstructorsData.get thy) rname)
-         handle Option => raise Match;
+         handle Option.Option => raise Match;
        val new =
            if #big_rec_name lcon_info = #big_rec_name rcon_info
                andalso not (null (#free_iffs lcon_info)) then