src/HOL/Bali/WellType.thy
changeset 13462 56610e2ba220
parent 13384 a34e38154413
child 13524 604d0f3622d6
--- a/src/HOL/Bali/WellType.thy	Tue Aug 06 11:20:47 2002 +0200
+++ b/src/HOL/Bali/WellType.thy	Tue Aug 06 11:22:05 2002 +0200
@@ -620,7 +620,7 @@
      _ $ (Const ("Pair", _) $ _ $ (Const ("Pair", _) $ _ $
        x))) $ _ )) = is_Inj x
 in
-  make_simproc name lhs pred (thm name)
+  cond_simproc name lhs pred (thm name)
 end
 
 val wt_expr_proc  = wt_fun "wt_expr_eq"  "In1l" "\<exists>T.  U=Inl T  \<and> E,dt\<Turnstile>t\<Colon>-T"