src/HOL/Wellfounded.thy
changeset 61943 7fba644ed827
parent 61799 4cf66f21b764
child 61952 546958347e05
--- a/src/HOL/Wellfounded.thy	Sun Dec 27 21:46:36 2015 +0100
+++ b/src/HOL/Wellfounded.thy	Sun Dec 27 22:07:17 2015 +0100
@@ -32,7 +32,7 @@
 text\<open>Restriction to domain @{term A} and range @{term B}.  If @{term r} is
     well-founded over their intersection, then @{term "wf r"}\<close>
 lemma wfI: 
- "[| r \<subseteq> A <*> B; 
+ "[| r \<subseteq> A \<times> B; 
      !!x P. [|\<forall>x. (\<forall>y. (y,x) : r --> P y) --> P x;  x : A; x : B |] ==> P x |]
   ==>  wf r"
   unfolding wf_def by blast